src/HOL/ex/Reflection_Examples.thy
changeset 66453 cc19f7ca2ed6
parent 61933 cf58b5b794b2
child 69597 ff784d5a5bfb
equal deleted inserted replaced
66452:450cefec7c11 66453:cc19f7ca2ed6
     3 *)
     3 *)
     4 
     4 
     5 section \<open>Examples for generic reflection and reification\<close>
     5 section \<open>Examples for generic reflection and reification\<close>
     6 
     6 
     7 theory Reflection_Examples
     7 theory Reflection_Examples
     8 imports Complex_Main "~~/src/HOL/Library/Reflection"
     8 imports Complex_Main "HOL-Library.Reflection"
     9 begin
     9 begin
    10 
    10 
    11 text \<open>This theory presents two methods: reify and reflection\<close>
    11 text \<open>This theory presents two methods: reify and reflection\<close>
    12 
    12 
    13 text \<open>
    13 text \<open>