src/FOL/ex/Locale_Test/Locale_Test1.thy
changeset 67740 b6ce18784872
parent 67450 b0ae74b86ef3
child 69054 ba8104f79d7b
equal deleted inserted replaced
67739:e512938b853c 67740:b6ce18784872
   521   x.lor_triv
   521   x.lor_triv
   522 
   522 
   523 
   523 
   524 subsection \<open>Rewrite morphisms in expressions\<close>
   524 subsection \<open>Rewrite morphisms in expressions\<close>
   525 
   525 
   526 interpretation y: logic_o "(\<or>)" "Not" replaces bool_logic_o2: "logic_o.lor_o((\<or>), Not, x, y) \<longleftrightarrow> x \<and> y"
   526 interpretation y: logic_o "(\<or>)" "Not" rewrites bool_logic_o2: "logic_o.lor_o((\<or>), Not, x, y) \<longleftrightarrow> x \<and> y"
   527 proof -
   527 proof -
   528   show bool_logic_o: "PROP logic_o((\<or>), Not)" by unfold_locales fast+
   528   show bool_logic_o: "PROP logic_o((\<or>), Not)" by unfold_locales fast+
   529   show "logic_o.lor_o((\<or>), Not, x, y) \<longleftrightarrow> x \<and> y" unfolding logic_o.lor_o_def [OF bool_logic_o] by fast
   529   show "logic_o.lor_o((\<or>), Not, x, y) \<longleftrightarrow> x \<and> y" unfolding logic_o.lor_o_def [OF bool_logic_o] by fast
   530 qed
   530 qed
   531 
   531