src/HOL/MicroJava/DFA/Semilattices.thy
author paulson <lp15@cam.ac.uk>
Wed, 01 Apr 2015 16:04:21 +0100
changeset 59872 db4000b71fdb
parent 58886 8a6cac7c7247
child 61361 8b5f00202e1a
permissions -rw-r--r--
Theorem "arctan" is no longer a default simprule

(*  Title:      HOL/MicroJava/DFA/Semilattices.thy
    Author:     Gerwin Klein
    Copyright   2003 TUM
*)

section {* Semilattices *}

(*<*)
theory Semilattices
imports Err Opt Product Listn
begin

end
(*>*)