src/FOL/ex/LocaleTest.thy
changeset 24788 f0dba1cda0b5
parent 24499 5a3ee202e0b0
child 25282 1cc04c8e1253
equal deleted inserted replaced
24787:df56433cc059 24788:f0dba1cda0b5
   207   print_interps! IA
   207   print_interps! IA
   208   fix beta and gamma
   208   fix beta and gamma
   209   interpret i9: ID [a beta _]
   209   interpret i9: ID [a beta _]
   210     apply - apply assumption
   210     apply - apply assumption
   211     apply unfold_locales
   211     apply unfold_locales
       
   212     apply (rule refl) (*FIXME: should have been discharged by unfold_locales*)
   212     apply (rule refl) done
   213     apply (rule refl) done
   213 qed rule
   214 qed rule
   214 
   215 
   215 
   216 
   216 (* Definition involving free variable *)
   217 (* Definition involving free variable *)