src/HOL/Finite_Set.thy
changeset 15770 90b6433c6093
parent 15765 6472d4942992
child 15780 6744bba5561d
equal deleted inserted replaced
15769:38c8ea8521e7 15770:90b6433c6093
  2306 using Distrib_Lattice_min_max
  2306 using Distrib_Lattice_min_max
  2307 by (fast dest: Distrib_Lattice.axioms)
  2307 by (fast dest: Distrib_Lattice.axioms)
  2308 
  2308 
  2309 text {* Classical rules from the locales are deleted in the above
  2309 text {* Classical rules from the locales are deleted in the above
  2310   interpretations, since they interfere with the claset setup for
  2310   interpretations, since they interfere with the claset setup for
  2311   {text "op \<le>"}. *)
  2311   @{text "op \<le>"}. *}
  2312 
  2312 
  2313 text{* Now we instantiate the recursion equations and declare them
  2313 text{* Now we instantiate the recursion equations and declare them
  2314 simplification rules: *}
  2314 simplification rules: *}
  2315 
  2315 
  2316 (* Making Min (resp. Max) a defined parameter of a locale suitably
  2316 (* Making Min (resp. Max) a defined parameter of a locale suitably