(* * Copyright 2016, NICTA * * This software may be distributed and modified according to the terms of * the BSD 2-Clause license. Note that NO WARRANTY is provided. * See "LICENSE_BSD2.txt" for details. * * @TAG(NICTA_BSD) *) theory ShowTypes_Test imports Lib.ShowTypes CLib.LemmaBucket_C CParser.CTranslation begin text \ Simple demo and test. The main HOL theories don't have that much hidden polymorphism, so we use l4.verified. \ experiment begin lemma c_guard_cast_byte: "c_guard (x :: ('a :: {mem_type}) ptr) \ c_guard (ptr_coerce x :: 8 word ptr)" goal_show_types 0 using [[show_sorts]] goal_show_types 0 apply (case_tac x) apply (fastforce intro!: byte_ptr_guarded simp: c_guard_def dest: c_null_guard) done thm c_guard_cast_byte[where x = "Ptr (ucast (0 :: 8 word))"] thm_show_types c_guard_cast_byte[where x = "Ptr (ucast (0 :: 8 word))"] (* Round-trip test *) ML \ let val ctxt = Config.put show_sorts true @{context} (* NB: this test fails if we leave some polymorphism in the term *) val term = @{thm c_guard_cast_byte[where x = "Ptr (ucast (0 :: 8 word)) :: unit ptr"]} |> Thm.prop_of val string_no_types = Syntax.pretty_term ctxt term |> Pretty.string_of |> YXML.content_of val string_show_types = Show_Types.term_show_types true ctxt term val _ = assert (Syntax.read_term ctxt string_no_types <> term) "Show_Types test (baseline)" val _ = assert (Syntax.read_term ctxt string_show_types = term) "Show_Types test" in () end \ end end